Skip to content
This repository has been archived by the owner on Sep 25, 2020. It is now read-only.

Protocol_Main breaks simplifier #61

Closed
dominique-unruh opened this issue Jul 9, 2017 · 2 comments
Closed

Protocol_Main breaks simplifier #61

dominique-unruh opened this issue Jul 9, 2017 · 2 comments

Comments

@dominique-unruh
Copy link
Contributor

In the following code, the by simp command fails, even though test_def is a simplifier rule.
When replacing imports Protocol_Main by imports Main, the by simp command works.
(This problem also occurs when one programatically access the simplifier via libisabelle.)

theory Scratch  
  imports Protocol_Main
begin
  
definition test where "test (x::int) = x"
declare test_def[simp]
  
lemma test2: "a=1 ⟶ test a=1"
  by simp 
@larsrh
Copy link
Owner

larsrh commented Jul 10, 2017

I vaguely remember this problem from updating Leon to Isabelle2016-1. The solution is to reorder imports in Protocol_Main. I'll try to fix this today and push out a new release.

@larsrh larsrh closed this as completed in eaafee2 Jul 10, 2017
@larsrh
Copy link
Owner

larsrh commented Jul 10, 2017

Fixed in 0.8.3.

Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
None yet
Projects
None yet
Development

No branches or pull requests

2 participants