src/HOL/Tools/Nitpick/nitpick_hol.ML
changeset 56245 84fc7dfa3cd4
parent 56243 2e10a36b8d46
child 57227 4c2156fdfe71
--- a/src/HOL/Tools/Nitpick/nitpick_hol.ML	Fri Mar 21 15:12:03 2014 +0100
+++ b/src/HOL/Tools/Nitpick/nitpick_hol.ML	Fri Mar 21 20:33:56 2014 +0100
@@ -363,9 +363,9 @@
    "Nitpick_Nut.nut_from_term", and perhaps in "Nitpick_Mono.consider_term" as
    well. *)
 val built_in_consts =
-  [(@{const_name all}, 1),
-   (@{const_name "=="}, 2),
-   (@{const_name "==>"}, 2),
+  [(@{const_name Pure.all}, 1),
+   (@{const_name Pure.eq}, 2),
+   (@{const_name Pure.imp}, 2),
    (@{const_name Pure.conjunction}, 2),
    (@{const_name Trueprop}, 1),
    (@{const_name Not}, 1),
@@ -973,7 +973,7 @@
       fold (fn (z as ((s, _), T)) => fn t' =>
                Logic.all_const T $ Abs (s, T, abstract_over (Var z, t')))
            (take (length zs' - length zs) zs')
-    fun aux zs (@{const "==>"} $ t1 $ t2) =
+    fun aux zs (@{const Pure.imp} $ t1 $ t2) =
         let val zs' = Term.add_vars t1 zs in
           close_up zs zs' (Logic.mk_implies (t1, aux zs' t2))
         end
@@ -1178,7 +1178,7 @@
   | loose_bvar1_count (Abs (_, _, t), k) = loose_bvar1_count (t, k + 1)
   | loose_bvar1_count _ = 0
 
-fun s_betapply _ (t1 as Const (@{const_name "=="}, _) $ t1', t2) =
+fun s_betapply _ (t1 as Const (@{const_name Pure.eq}, _) $ t1', t2) =
     if t1' aconv t2 then @{prop True} else t1 $ t2
   | s_betapply _ (t1 as Const (@{const_name HOL.eq}, _) $ t1', t2) =
     if t1' aconv t2 then @{term True} else t1 $ t2
@@ -1422,8 +1422,8 @@
    simplification rules (equational specifications). *)
 fun term_under_def t =
   case t of
-    @{const "==>"} $ _ $ t2 => term_under_def t2
-  | Const (@{const_name "=="}, _) $ t1 $ _ => term_under_def t1
+    @{const Pure.imp} $ _ $ t2 => term_under_def t2
+  | Const (@{const_name Pure.eq}, _) $ t1 $ _ => term_under_def t1
   | @{const Trueprop} $ t1 => term_under_def t1
   | Const (@{const_name HOL.eq}, _) $ t1 $ _ => term_under_def t1
   | Abs (_, _, t') => term_under_def t'
@@ -1448,7 +1448,7 @@
       | aux _ _ = NONE
     val (lhs, rhs) =
       case t of
-        Const (@{const_name "=="}, _) $ t1 $ t2 => (t1, t2)
+        Const (@{const_name Pure.eq}, _) $ t1 $ t2 => (t1, t2)
       | @{const Trueprop} $ (Const (@{const_name HOL.eq}, _) $ t1 $ t2) =>
         (t1, t2)
       | _ => raise TERM ("Nitpick_HOL.normalized_rhs_of", [t])
@@ -1527,9 +1527,9 @@
 
 fun lhs_of_equation t =
   case t of
-    Const (@{const_name all}, _) $ Abs (_, _, t1) => lhs_of_equation t1
-  | Const (@{const_name "=="}, _) $ t1 $ _ => SOME t1
-  | @{const "==>"} $ _ $ t2 => lhs_of_equation t2
+    Const (@{const_name Pure.all}, _) $ Abs (_, _, t1) => lhs_of_equation t1
+  | Const (@{const_name Pure.eq}, _) $ t1 $ _ => SOME t1
+  | @{const Pure.imp} $ _ $ t2 => lhs_of_equation t2
   | @{const Trueprop} $ t1 => lhs_of_equation t1
   | Const (@{const_name All}, _) $ Abs (_, _, t1) => lhs_of_equation t1
   | Const (@{const_name HOL.eq}, _) $ t1 $ _ => SOME t1
@@ -1947,7 +1947,7 @@
           @{const Trueprop} $ extensional_equal j T t1 t2
         | @{const Trueprop} $ t' =>
           @{const Trueprop} $ HOLogic.mk_eq (t', @{const True})
-        | Const (@{const_name "=="}, Type (_, [T, _])) $ t1 $ t2 =>
+        | Const (@{const_name Pure.eq}, Type (_, [T, _])) $ t1 $ t2 =>
           @{const Trueprop} $ extensional_equal j T t1 t2
         | _ => (warning ("Ignoring " ^ quote tag ^ " for non-equation " ^
                          quote (Syntax.string_of_term ctxt t) ^ ".");