src/HOL/Decision_Procs/Commutative_Ring.thy
changeset 47432 e1576d13e933
parent 41807 ab5d2d81f9fb
child 48891 c0eafbd55de3
equal deleted inserted replaced
47431:d9dd4a9f18fc 47432:e1576d13e933
   312   then show ?thesis by (simp only: norm_ci)
   312   then show ?thesis by (simp only: norm_ci)
   313 qed
   313 qed
   314 
   314 
   315 
   315 
   316 use "commutative_ring_tac.ML"
   316 use "commutative_ring_tac.ML"
   317 setup Commutative_Ring_Tac.setup
   317 
       
   318 method_setup comm_ring = {*
       
   319   Scan.succeed (SIMPLE_METHOD' o Commutative_Ring_Tac.tac)
       
   320 *} "reflective decision procedure for equalities over commutative rings"
   318 
   321 
   319 end
   322 end