src/HOL/ex/MT.thy
changeset 3842 b55686a7b22c
parent 1476 608483c2122a
child 5102 8c782c25a11e
--- a/src/HOL/ex/MT.thy	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOL/ex/MT.thy	Fri Oct 10 19:02:28 1997 +0200
@@ -247,7 +247,7 @@
      ve_dom(ve) = te_dom(te) & 
      ( ! x. 
          x:ve_dom(ve) --> 
-         (? c.ve_app ve x = v_const(c) & c isof te_app te x) 
+         (? c. ve_app ve x = v_const(c) & c isof te_app te x) 
      ) 
    "
 
@@ -263,7 +263,7 @@
            p = (v_clos(<|ev,e,ve|>),t) & 
            te |- fn ev => e ===> t & 
            ve_dom(ve) = te_dom(te) & 
-           (! ev1.ev1:ve_dom(ve) --> (ve_app ve ev1,te_app te ev1) : r) 
+           (! ev1. ev1:ve_dom(ve) --> (ve_app ve ev1,te_app te ev1) : r) 
        ) 
      } 
    "