src/HOL/HOL.thy
changeset 22993 838c66e760b5
parent 22839 ede26eb5e549
child 23037 6c72943a71b1
--- a/src/HOL/HOL.thy	Thu May 17 19:29:39 2007 +0200
+++ b/src/HOL/HOL.thy	Thu May 17 19:49:16 2007 +0200
@@ -227,7 +227,7 @@
   fun tr' c = (c, fn show_sorts => fn T => fn ts =>
     if T = dummyT orelse not (! show_types) andalso can Term.dest_Type T then raise Match
     else Syntax.const Syntax.constrainC $ Syntax.const c $ Syntax.term_of_typ show_sorts T);
-in map tr' [@{const_syntax "HOL.one"}, @{const_syntax "HOL.zero"}] end;
+in map tr' [@{const_syntax HOL.one}, @{const_syntax HOL.zero}] end;
 *} -- {* show types that are presumably too general *}
 
 
@@ -913,7 +913,7 @@
 struct
   type claset = Classical.claset
   val equality_name = @{const_name "op ="}
-  val not_name = @{const_name "Not"}
+  val not_name = @{const_name Not}
   val notE = @{thm HOL.notE}
   val ccontr = @{thm HOL.ccontr}
   val contr_tac = Classical.contr_tac