]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/assembly/compiler/tests.ma
mod change (-x)
[helm.git] / helm / software / matita / contribs / assembly / compiler / tests.ma
old mode 100755 (executable)
new mode 100644 (file)
index e07e440..344ac7c
@@ -225,4 +225,5 @@ lemma pippo : ∃b.preast_to_ast parsingResult = Some ? b.
  exists;
  [ apply (match preast_to_ast parsingResult with [ None ⇒ AST_ROOT (AST_NO_DECL O empty_env []) | Some x ⇒ x]);
  | reflexivity
- ].
+ ]
+qed.