schematic goals;
authorwenzelm
Fri, 01 Dec 2000 19:42:05 +0100
changeset 10567 e7c9900cca4d
parent 10566 7ed4f5a6c63f
child 10568 a7701b1d6c6a
schematic goals;
src/HOL/Lambda/Type.thy
--- a/src/HOL/Lambda/Type.thy	Fri Dec 01 19:41:45 2000 +0100
+++ b/src/HOL/Lambda/Type.thy	Fri Dec 01 19:42:05 2000 +0100
@@ -59,16 +59,12 @@
 
 subsection {* Some examples *}
 
-lemma "\<exists>T U. e |- Abs (Abs (Abs (Var 1 $ (Var 2 $ Var 1 $ Var 0)))) : T \<and> U = T"
-  apply (intro exI conjI)
-   apply force
-  apply (rule refl)
+lemma "e |- Abs (Abs (Abs (Var 1 $ (Var 2 $ Var 1 $ Var 0)))) : ?T"
+  apply force
   done
 
-lemma "\<exists>T U. e |- Abs (Abs (Abs (Var 2 $ Var 0 $ (Var 1 $ Var 0)))) : T \<and> U = T";
-  apply (intro exI conjI)
-   apply force
-  apply (rule refl)
+lemma "e |- Abs (Abs (Abs (Var 2 $ Var 0 $ (Var 1 $ Var 0)))) : ?T"
+  apply force
   done